aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/Sendback.thy
blob: f14ae72c2530e3293c410abb3f6997aef26d22e6 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
(* Demonstrate the use of literal command markup *)

theory Sendback imports Main begin

ML {* val pgasciiN = "PGASCII";
fun special oct =
  if print_mode_active pgasciiN then chr 1 ^ chr (ord (oct_char oct) - 167)
  else oct_char oct; 
fun sendback cmd = writeln ("Try this: \n   " ^ (special "375") ^ cmd ^ "\n\n")
*}

theorem and_comms: "A & B --> B & A"
proof
  ML {* sendback "assume \"A & B\"" *}
  ML {* sendback "then; show \"B & A\"" *}
  ML {* sendback "proof; assume B and A; then" *}
  ML {* sendback "show ?thesis; ..; qed" *}
  ML {* sendback "qed" *}
qed