--- a/src/CCL/CCL.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/CCL/CCL.thy Wed Apr 28 12:07:52 2010 +0200
@@ -17,7 +17,7 @@
*}
classes prog < "term"
-defaultsort prog
+default_sort prog
arities "fun" :: (prog, prog) prog
--- a/src/FOL/IFOL.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/FOL/IFOL.thy Wed Apr 28 12:07:52 2010 +0200
@@ -31,7 +31,7 @@
global
classes "term"
-defaultsort "term"
+default_sort "term"
typedecl o
--- a/src/FOLP/IFOLP.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/FOLP/IFOLP.thy Wed Apr 28 12:07:52 2010 +0200
@@ -15,7 +15,7 @@
global
classes "term"
-defaultsort "term"
+default_sort "term"
typedecl p
typedecl o
--- a/src/HOL/HOL.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOL/HOL.thy Wed Apr 28 12:07:52 2010 +0200
@@ -40,7 +40,7 @@
subsubsection {* Core syntax *}
classes type
-defaultsort type
+default_sort type
setup {* Object_Logic.add_base_sort @{sort type} *}
arities
--- a/src/HOL/ex/Higher_Order_Logic.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOL/ex/Higher_Order_Logic.thy Wed Apr 28 12:07:52 2010 +0200
@@ -20,7 +20,7 @@
subsection {* Pure Logic *}
classes type
-defaultsort type
+default_sort type
typedecl o
arities
--- a/src/HOLCF/Adm.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Adm.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Cont
begin
-defaultsort cpo
+default_sort cpo
subsection {* Definitions *}
--- a/src/HOLCF/Algebraic.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Algebraic.thy Wed Apr 28 12:07:52 2010 +0200
@@ -297,7 +297,7 @@
subsection {* Type constructor for finite deflations *}
-defaultsort profinite
+default_sort profinite
typedef (open) 'a fin_defl = "{d::'a \<rightarrow> 'a. finite_deflation d}"
by (fast intro: finite_deflation_approx)
--- a/src/HOLCF/Cfun.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Cfun.thy Wed Apr 28 12:07:52 2010 +0200
@@ -9,7 +9,7 @@
imports Pcpodef Ffun Product_Cpo
begin
-defaultsort cpo
+default_sort cpo
subsection {* Definition of continuous function type *}
@@ -511,7 +511,7 @@
subsection {* Strictified functions *}
-defaultsort pcpo
+default_sort pcpo
definition
strictify :: "('a \<rightarrow> 'b) \<rightarrow> 'a \<rightarrow> 'b" where
--- a/src/HOLCF/CompactBasis.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/CompactBasis.thy Wed Apr 28 12:07:52 2010 +0200
@@ -10,7 +10,7 @@
subsection {* Compact bases of bifinite domains *}
-defaultsort profinite
+default_sort profinite
typedef (open) 'a compact_basis = "{x::'a::profinite. compact x}"
by (fast intro: compact_approx)
--- a/src/HOLCF/Cont.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Cont.thy Wed Apr 28 12:07:52 2010 +0200
@@ -14,7 +14,7 @@
of default class po
*}
-defaultsort po
+default_sort po
subsection {* Definitions *}
--- a/src/HOLCF/Cprod.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Cprod.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Bifinite
begin
-defaultsort cpo
+default_sort cpo
subsection {* Continuous case function for unit type *}
--- a/src/HOLCF/Deflation.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Deflation.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Cfun
begin
-defaultsort cpo
+default_sort cpo
subsection {* Continuous deflations *}
--- a/src/HOLCF/Domain.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Domain.thy Wed Apr 28 12:07:52 2010 +0200
@@ -16,7 +16,7 @@
("Tools/Domain/domain_extender.ML")
begin
-defaultsort pcpo
+default_sort pcpo
subsection {* Casedist *}
--- a/src/HOLCF/FOCUS/Fstream.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/FOCUS/Fstream.thy Wed Apr 28 12:07:52 2010 +0200
@@ -12,7 +12,7 @@
imports "../ex/Stream"
begin
-defaultsort type
+default_sort type
types 'a fstream = "'a lift stream"
--- a/src/HOLCF/FOCUS/Fstreams.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/FOCUS/Fstreams.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
theory Fstreams imports "../ex/Stream" begin
-defaultsort type
+default_sort type
types 'a fstream = "('a lift) stream"
--- a/src/HOLCF/Fix.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Fix.thy Wed Apr 28 12:07:52 2010 +0200
@@ -9,7 +9,7 @@
imports Cfun
begin
-defaultsort pcpo
+default_sort pcpo
subsection {* Iteration *}
--- a/src/HOLCF/Fixrec.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Fixrec.thy Wed Apr 28 12:07:52 2010 +0200
@@ -13,7 +13,7 @@
subsection {* Maybe monad type *}
-defaultsort cpo
+default_sort cpo
pcpodef (open) 'a maybe = "UNIV::(one ++ 'a u) set"
by simp_all
@@ -463,7 +463,7 @@
subsection {* Match functions for built-in types *}
-defaultsort pcpo
+default_sort pcpo
definition
match_UU :: "'a \<rightarrow> 'c maybe \<rightarrow> 'c maybe"
--- a/src/HOLCF/HOLCF.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/HOLCF.thy Wed Apr 28 12:07:52 2010 +0200
@@ -12,7 +12,7 @@
Sum_Cpo
begin
-defaultsort pcpo
+default_sort pcpo
text {* Legacy theorem names *}
--- a/src/HOLCF/IOA/Storage/Correctness.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/Storage/Correctness.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports SimCorrectness Spec Impl
begin
-defaultsort type
+default_sort type
definition
sim_relation :: "((nat * bool) * (nat set * bool)) set" where
--- a/src/HOLCF/IOA/meta_theory/Abstraction.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Abstraction.thy Wed Apr 28 12:07:52 2010 +0200
@@ -9,7 +9,7 @@
uses ("automaton.ML")
begin
-defaultsort type
+default_sort type
definition
cex_abs :: "('s1 => 's2) => ('a,'s1)execution => ('a,'s2)execution" where
--- a/src/HOLCF/IOA/meta_theory/Automata.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Automata.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Asig
begin
-defaultsort type
+default_sort type
types
('a, 's) transition = "'s * 'a * 's"
--- a/src/HOLCF/IOA/meta_theory/LiveIOA.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/LiveIOA.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports TLS
begin
-defaultsort type
+default_sort type
types
('a, 's) live_ioa = "('a,'s)ioa * ('a,'s)ioa_temp"
--- a/src/HOLCF/IOA/meta_theory/Pred.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Pred.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Main
begin
-defaultsort type
+default_sort type
types
'a predicate = "'a => bool"
--- a/src/HOLCF/IOA/meta_theory/RefMappings.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/RefMappings.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Traces
begin
-defaultsort type
+default_sort type
definition
move :: "[('a,'s)ioa,('a,'s)pairs,'s,'a,'s] => bool" where
--- a/src/HOLCF/IOA/meta_theory/Sequence.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Sequence.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Seq
begin
-defaultsort type
+default_sort type
types 'a Seq = "'a::type lift seq"
--- a/src/HOLCF/IOA/meta_theory/Simulations.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Simulations.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports RefCorrectness
begin
-defaultsort type
+default_sort type
definition
is_simulation :: "[('s1 * 's2)set,('a,'s1)ioa,('a,'s2)ioa] => bool" where
--- a/src/HOLCF/IOA/meta_theory/TL.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/TL.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Pred Sequence
begin
-defaultsort type
+default_sort type
types
'a temporal = "'a Seq predicate"
--- a/src/HOLCF/IOA/meta_theory/TLS.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/TLS.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports IOA TL
begin
-defaultsort type
+default_sort type
types
('a, 's) ioa_temp = "('a option,'s)transition temporal"
--- a/src/HOLCF/IOA/meta_theory/Traces.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Traces.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Sequence Automata
begin
-defaultsort type
+default_sort type
types
('a,'s)pairs = "('a * 's) Seq"
--- a/src/HOLCF/Lift.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Lift.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Discrete Up Countable
begin
-defaultsort type
+default_sort type
pcpodef 'a lift = "UNIV :: 'a discr u set"
by simp_all
--- a/src/HOLCF/Product_Cpo.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Product_Cpo.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Adm
begin
-defaultsort cpo
+default_sort cpo
subsection {* Unit type is a pcpo *}
--- a/src/HOLCF/Representable.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Representable.thy Wed Apr 28 12:07:52 2010 +0200
@@ -42,7 +42,7 @@
@{term rep}, unless specified otherwise.
*}
-defaultsort rep
+default_sort rep
subsection {* Representations of types *}
--- a/src/HOLCF/Sprod.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Sprod.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Bifinite
begin
-defaultsort pcpo
+default_sort pcpo
subsection {* Definition of strict product type *}
--- a/src/HOLCF/Ssum.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Ssum.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Tr
begin
-defaultsort pcpo
+default_sort pcpo
subsection {* Definition of strict sum type *}
--- a/src/HOLCF/Tr.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Tr.thy Wed Apr 28 12:07:52 2010 +0200
@@ -62,7 +62,7 @@
subsection {* Case analysis *}
-defaultsort pcpo
+default_sort pcpo
definition
trifte :: "'c \<rightarrow> 'c \<rightarrow> tr \<rightarrow> 'c" where
--- a/src/HOLCF/Universal.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Universal.thy Wed Apr 28 12:07:52 2010 +0200
@@ -340,7 +340,7 @@
subsection {* Universality of \emph{udom} *}
-defaultsort bifinite
+default_sort bifinite
subsubsection {* Choosing a maximal element from a finite set *}
--- a/src/HOLCF/Up.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/Up.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports Bifinite
begin
-defaultsort cpo
+default_sort cpo
subsection {* Definition of new type for lifting *}
--- a/src/HOLCF/ex/Domain_Proofs.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/ex/Domain_Proofs.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports HOLCF
begin
-defaultsort rep
+default_sort rep
(*
--- a/src/HOLCF/ex/Letrec.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/ex/Letrec.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports HOLCF
begin
-defaultsort pcpo
+default_sort pcpo
definition
CLetrec :: "('a \<rightarrow> 'a \<times> 'b) \<rightarrow> 'b" where
--- a/src/HOLCF/ex/New_Domain.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/ex/New_Domain.thy Wed Apr 28 12:07:52 2010 +0200
@@ -13,7 +13,7 @@
i.e. types in class @{text rep}.
*}
-defaultsort rep
+default_sort rep
text {*
Provided that @{text rep} is the default sort, the @{text new_domain}
--- a/src/HOLCF/ex/Powerdomain_ex.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/ex/Powerdomain_ex.thy Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
imports HOLCF
begin
-defaultsort bifinite
+default_sort bifinite
subsection {* Monadic sorting example *}
--- a/src/LCF/LCF.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/LCF/LCF.thy Wed Apr 28 12:07:52 2010 +0200
@@ -14,7 +14,7 @@
subsection {* Natural Deduction Rules for LCF *}
classes cpo < "term"
-defaultsort cpo
+default_sort cpo
typedecl tr
typedecl void
--- a/src/Pure/Isar/isar_syn.ML Wed Apr 28 11:41:27 2010 +0200
+++ b/src/Pure/Isar/isar_syn.ML Wed Apr 28 12:07:52 2010 +0200
@@ -96,7 +96,7 @@
>> (Toplevel.theory o AxClass.axiomatize_classrel_cmd));
val _ =
- OuterSyntax.local_theory "defaultsort" "declare default sort for explicit type variables"
+ OuterSyntax.local_theory "default_sort" "declare default sort for explicit type variables"
K.thy_decl
(P.sort >> (fn s => fn lthy => Local_Theory.set_defsort (Syntax.read_sort lthy s) lthy));
--- a/src/Sequents/LK0.thy Wed Apr 28 11:41:27 2010 +0200
+++ b/src/Sequents/LK0.thy Wed Apr 28 12:07:52 2010 +0200
@@ -15,7 +15,7 @@
global
classes "term"
-defaultsort "term"
+default_sort "term"
consts