aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/trac/trac-307.thy
blob: b4d69be23c356fd7064d3423e848946ce6cd205e (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15

theory trac307 imports Main begin

lemma foo: "Suc x = Suc x" ..

(* 2. Go to the simp-command that does not terminate
   3. Perform the following actions:
      Undo, Interrupt, Undo, Next
   Sync is lost.
*)

lemma "P (Suc x)" apply (simp add: foo)

end