diff -r 143f58bb34f9 -r 0909deb8059b src/HOL/Nominal/Examples/SOS.thy --- a/src/HOL/Nominal/Examples/SOS.thy Thu May 26 16:57:14 2016 +0200 +++ b/src/HOL/Nominal/Examples/SOS.thy Thu May 26 17:51:22 2016 +0200 @@ -16,7 +16,7 @@ atom_decl name -text {* types and terms *} +text \types and terms\ nominal_datatype ty = TVar "nat" | Arrow "ty" "ty" ("_\_" [100,100] 100) @@ -33,7 +33,7 @@ by (induct T rule: ty.induct) (auto simp add: fresh_nat) -text {* Parallel and single substitution. *} +text \Parallel and single substitution.\ fun lookup :: "(name\trm) list \ name \ trm" where @@ -94,7 +94,7 @@ by (nominal_induct t rule: trm.strong_induct) (auto simp add: fresh_list_nil) -text {* Single substitution *} +text \Single substitution\ abbreviation subst :: "trm \ name \ trm \ trm" ("_[_::=_]" [100,100,100] 100) where @@ -126,7 +126,7 @@ by (nominal_induct e avoiding: \ x e' rule: trm.strong_induct) (auto simp add: fresh_list_cons fresh_atm forget lookup_fresh lookup_fresh') -text {* Typing Judgements *} +text \Typing Judgements\ inductive valid :: "(name\ty) list \ bool" @@ -158,7 +158,7 @@ using a1 a2 a3 by (induct) (auto simp add: fresh_set fresh_prod fresh_atm) -text {* Typing Relation *} +text \Typing Relation\ inductive typing :: "(name\ty) list\trm\ty\bool" ("_ \ _ : _" [60,60,60] 60) @@ -244,7 +244,7 @@ using a b type_substitutivity_aux[where \="[]"] by (auto) -text {* Values *} +text \Values\ inductive val :: "trm\bool" where @@ -258,7 +258,7 @@ "\ val (Var x)" by (auto elim: val.cases) -text {* Big-Step Evaluation *} +text \Big-Step Evaluation\ inductive big :: "trm\trm\bool" ("_ \ _" [80,80] 80) @@ -428,7 +428,7 @@ shows "v \ v" using a by (simp add: values_reduce_to_themselves Vs_are_values) -text {* '\ maps x to e' asserts that \ substitutes x with e *} +text \'\ maps x to e' asserts that \ substitutes x with e\ abbreviation mapsto :: "(name\trm) list \ name \ trm \ bool" ("_ maps _ to _" [55,55,55] 55) where