src/HOL/Predicate.thy
changeset 23389 aaca6a8e5414
parent 22846 fb79144af9a3
child 23708 b5eb0b4dd17d
--- a/src/HOL/Predicate.thy	Thu Jun 14 18:33:29 2007 +0200
+++ b/src/HOL/Predicate.thy	Thu Jun 14 18:33:31 2007 +0200
@@ -34,11 +34,11 @@
 proof
   fix S
   assume "!!S. PROP P S"
-  show "PROP P (Collect S)" .
+  then show "PROP P (Collect S)" .
 next
   fix S
   assume "!!S. PROP P (Collect S)"
-  have "PROP P {x. x : S}" .
+  then have "PROP P {x. x : S}" .
   thus "PROP P S" by simp
 qed
 
@@ -46,11 +46,11 @@
 proof
   fix S
   assume "!!S. PROP P S"
-  show "PROP P (member S)" .
+  then show "PROP P (member S)" .
 next
   fix S
   assume "!!S. PROP P (member S)"
-  have "PROP P (member {x. S x})" .
+  then have "PROP P (member {x. S x})" .
   thus "PROP P S" by simp
 qed
 
@@ -96,11 +96,11 @@
 proof
   fix S
   assume "!!S. PROP P S"
-  show "PROP P (Collect2 S)" .
+  then show "PROP P (Collect2 S)" .
 next
   fix S
   assume "!!S. PROP P (Collect2 S)"
-  have "PROP P (Collect2 (member2 S))" .
+  then have "PROP P (Collect2 (member2 S))" .
   thus "PROP P S" by simp
 qed
 
@@ -108,11 +108,11 @@
 proof
   fix S
   assume "!!S. PROP P S"
-  show "PROP P (member2 S)" .
+  then show "PROP P (member2 S)" .
 next
   fix S
   assume "!!S. PROP P (member2 S)"
-  have "PROP P (member2 (Collect2 S))" .
+  then have "PROP P (member2 (Collect2 S))" .
   thus "PROP P S" by simp
 qed