src/HOLCF/IOA/NTP/Lemmas.ML
changeset 4423 a129b817b58a
parent 4377 2cba48b0f1c4
child 4532 006e5572aca8
--- a/src/HOLCF/IOA/NTP/Lemmas.ML	Tue Dec 16 15:17:26 1997 +0100
+++ b/src/HOLCF/IOA/NTP/Lemmas.ML	Tue Dec 16 17:58:03 1997 +0100
@@ -7,7 +7,7 @@
 
 (* Logic *)
 val prems = goal HOL.thy "(P ==> Q-->R) ==> P&Q --> R";
-  by(fast_tac (claset() addDs prems) 1);
+  by (fast_tac (claset() addDs prems) 1);
 qed "imp_conj_lemma";
 
 goal HOL.thy "(A --> B & C) = ((A --> B) & (A --> C))";
@@ -35,8 +35,8 @@
 (* Arithmetic *)
 
 goal Arith.thy "!!x. 0<x ==> (x-1 = y) = (x = Suc(y))";
-by(asm_simp_tac (simpset() addsimps [diff_Suc] addsplits [expand_nat_case]) 1);
-by(Blast_tac 1);
+by (asm_simp_tac (simpset() addsimps [diff_Suc] addsplits [expand_nat_case]) 1);
+by (Blast_tac 1);
 qed "pred_suc";