Coq/SSReflect/MathComp による定理証明 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

Size: px
Start display at page:

Download "Coq/SSReflect/MathComp による定理証明 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです."

Transcription

1

2 Coq/SSReflect/MathComp による定理証明 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

3

4 i Coq/SS- Reflect/MathComp 1 1 Coq/SSReflect/MathComp

5 ii 1 Coq/SSReflect/MathComp

6 iii 1 Coq/SSReflect/MathComp Coq/SSReflect/MathComp Microsoft Windows Coq/SSReflect/MathComp move=>, move:, move: =>, move/ apply, apply=>, apply:, apply: =>, apply/ case, case:, case=>, case: =>, case=> [ ], case/ elim, elim:, elim=>, elim: =>, elim=> [ ] rewrite move/, apply/, case/ have suff wlog Definition, Lemma, Theorem, Corollary, Fact, Proposition, Remark, Proof, Qed, Fixpoint Compute Check About Print Search Locate Abort Admitted Variable(s) Hypothesis Axiom Inductive 117

7 iv 3.15 Record Canonical Coq split left right exists MathComp ssrbool.v bool eqtype.v eqtype ssrnat.v SSReflect nat seq.v seq fintype.v bigop.v fintype finset Infotheo

8 1 1 Coq/SSReflect/MathComp Coq SSReflect MathComp Coq/SSReflect/MathComp

9 2 1 Coq/SSReflect/MathComp 1.1 Coq/SSReflect 1 /MathComp 1 Coq SSReflect MathComp Coq/SSReflect/ MathComp Coq/SSReflect/MathComp Coq/SSReflect/MathComp SSReflect 2 SSReflect Coq 1.1 Coq move=> A B C. forall A B C : Prop, (A -> B) /\ (B -> C) -> (A -> C) move=> A B C. A, B, C : Prop (A -> B) /\ (B -> C) -> (A -> C) 1.1 move=> A B C 1 2 Ssreflect Small Scale Reflection SSReflect

10 SSReflect A, B, C (A B) (B C) (A C) SSReflect forall A B C : Prop, (A -> B) /\ (B -> C) -> (A -> C). Proof. A, B, C move=> A B C. (A B) (B C) (A B) (B C) A B Hyp1 B C Hyp2 A C A Hyp3 C Hyp2 B B Hyp1 A A Hyp3 case. move=> Hyp1. move=> Hyp2. move=> Hyp3. apply: Hyp2. apply: Hyp1. by []. Qed. SSReflect 1.1 SSReflect SSReflect

11 4 1 Coq/SSReflect/MathComp Coq SSReflect INRIA Coq/SSReflect 15 7 MathComp Coq SSReflect 2 Coq, SSReflect Coq ACM (Association for Computing Machinery) 2013 ACM ACM SIGPLAN SSReflect 2011 EADS Georges Gonthier, 1962 Vladimir Voevodsky, EADS

12 Flyspeck Formal Proof of Kepler Conjecture IT C CompCert sel4 1 2 Johannes Kepler, Thomas Hales, 1958

13 6 1 Coq/SSReflect/MathComp Coq/SSReflect/MathComp ICT

14 1.2 7 Coq/SSReflect Coq/SSReflect Coq Coq Mizar 1 HOL Light 2 Agda Isabelle 3 Mizar a : A A a Mizar: HOL Light: Isabelle: Ernst Zermelo, Bertrand Russell, int, float

15 8 1 Coq/SSReflect/MathComp a A a A a A 1 a : A A a A B 1.2 A B A + B A B A B Σx : A, B A B A B Πx : A, B A B x A, B(x) Πx : A, B(x) A x B(x) x A, B(x) Σx : A, B(x) A x B(x) A B A + B A + B A B A + B A B A + B A B A B A + B B + A B + A b : B a : A A B Σx : A, B Σx : A, B (a, b) a : A b : B A B A, B A B A, B Σx : A, B Σx : A, B A, B A B 1 a A a : A a i A int i : int

16 25 2 Coq/SSReflect/MathComp Coq/SSReflect/MathComp

17 Coq 2.1 CoqIDE Proof General Coq Coq 2.1 P, Q : Prop Hyp : P P Q Prop Hyp P -> forall 1 -> 2.1 (P -> Q) -> P (P -> Q), P 2.1 1

18 Coq/SSReflect/MathComp Coq/SSReflect/MathComp CoqIDE From mathcomp Require Import ssreflect. Section ModusPonens. Variables X Y : Prop. Hypothesis XtoY_is_true : X -> Y. Hypothesis X_is_true : X. Theorem MP : Y. Proof. move: X_is_true. by []. Qed. End ModusPonens. Coq CoqIDE Coq 1 Coq 1

19 CoqIDE [Loading ML file ssreflect.cmxs... done] Coq SSReflect From mathcomp Require Import mathcomp ssreflect Coq SSReflect ssreflect div From mathcomp Require Import ssreflect div. From mathcomp Require Import ssreflect. From mathcomp Require Import div. 1 Section ModusPonens. Section ModusPonens End 1 Variables X Y : Prop. X is assumed Y is assumed

20 Variables 1 ModusPonens X, Y Variable Variable :. Variables... :. 2 X Y Prop Coq/SSReflect/MathComp 1 Hypothesis XtoY_is_true : X -> Y. XtoY_is_true is assumed Hypothesis X -> Y XtoY_is_true X Y > -> - > Coq X -> Y X -> Y X -> Y 1 X X_is_true 1 Theorem MP : Y. 1 2 Variables Variable Coq Variable Variables A E Variables A B... E Variables A B C D E

21 subgoal X, Y : Prop XtoY_is_true : X -> Y X_is_true : X (1/1) Y 1 Theorem Theorem... :. MP Y subgoal Theorem 4 subgoals X, Y : Prop X Y Prop Variable XtoY_is_true : X -> Y X_is_true : X Hypothesis (1/1) n / m 2.1 Coq X, Y : Prop XtoY_is_true : X -> Y X_is_true : X Y X, Y X Y X Y 1 Coq

22 SSReflect

23 From mathcomp 2 Require Import all_ssreflect. 3 4 Set Implicit Arguments. 5 Unset Strict Implicit. 6 Import Prenex Implicits. 1 2 MathComp SSReflect Coq 7 8 Definition myset (M : Type) := M -> Prop. 9 Definition belong {M : Type} (A : myset M) (x : M) : 10 Prop := A x. 11 Notation "x A" := (belong A x) (at level 11). 12 Axiom axiom_myset : forall (M : Type )( A : myset M), 13 forall (x : M), (x A) \/ ~(x A). x Coq/SSReflect M : Type mother set M M M -> Prop myset M myset M M -> Prop Coq Coq Sets.Ensembles Ensemble M A : myset M

24 x : M A A x (A x) belong A x A x : Prop x A belong A x A x : Prop belong { } {M : Type} { } Coq myset (M : Type) := M -> Prop x x A x / A myset T axiom_myset Definition myemptyset {M : Type} : myset M := fun _ => False. 16 Definition mymotherset {M : Type} : myset M := fun _ => True. myemptyset mymotherset x : M (x myemptyset) x : M x mymotherset 5.2 A, B A B x A x B mysub M -> mysub M -> Prop mysub M Prop mysub Definition mysub {M} := fun (A B : myset M) => 19 (forall (x : M), (x A) -> (x B)). 20 Notation "A B" := (mysub A B) (at level 11).

25 Section. 23 Variable M : Type Lemma Sub_Mother (A : myset M) : A mymotherset. 26 Proof. by []. Qed Lemma Sub_Empty (A : myset M) : myemptyset A. 29 Proof. by []. Qed Lemma rfl_sub (A : myset M) : (A A). 32 Proof. by []. Qed Lemma transitive_sub (A B C : myset M): 35 (A B) -> (B C) -> (A C). 36 Proof. by move=> H1 H2 t H3; apply: H2; apply: H1. Qed End. 2 Section M : Type Variable mysub Sub Sub_Mother mysub mymotherset Sub_Empty rfl_sub reflexivity rfl transitive_sub 1 A, B A = B A B B A Coq myset {M : Type} A = B A B B A

26 rewrite rfl_sub Definition eqmyset {M : Type }:= 41 fun (A B : myset M) => (A B /\ B A). 42 Axiom axiom_exteqmyset : forall {M : Type} (A B : myset M), 43 eqmyset A B -> A = B. axiom_exteqmyset Section. 46 Variable Mother : Type Lemma rfl_eqs (A : myset Mother) : A = A. 49 Proof. by []. Qed Lemma sym_eqs (A B : myset Mother) : A = B -> B = A. 52 Proof. move=> H. by rewrite H. Qed End. eq S myset eqs sym symmetry Definition mycomplement {M : Type} (A : myset M) : myset M := 57 fun (x : M) => ~(A x). 58 Notation "A ^c" := ( mycomplement A) (at level 11) Definition mycup {M : Type} (A B : myset M) : myset M := 61 fun (x : M) => (x A) \/ (x B). 62 Notation "A B" := (mycup A B) (at level 11). mycomplement A x A c

27 162 5 mycup \/ A B Section. 65 Variable M : Type Lemma cempty_mother : (@myemptyset M)^c = mymotherset. 68 Proof. 69 apply: axiom_exteqmyset; rewrite / eqmyset. 70 by apply: conj; rewrite / mysub / mycomplement // => x Hfull. 71 Qed Lemma cc_cancel (A : myset M) : (A^c)^c = A. 74 apply: axiom_exteqmyset; rewrite / eqmyset. 75 apply: conj; rewrite / mysub / mycomplement => x H //. 76 by case: ( axiom_myset A x). 77 Qed Lemma cmother_empty : (@mymotherset M)^c = myemptyset. 80 Proof. by rewrite - cempty_mother cc_cancel. Qed. M Coq Error: Cannot infer the implicit parameter M of mycomplement whose type is "Type" in environment: M : Type M myemptyset M M M Coq Lemma mycupa (A B C : myset M) : (A B) C = A (B C). 83 Proof.

28 apply: axiom_exteqmyset. 85 rewrite / eqmyset / mysub. 86 apply: conj => x [H1 H2]. 87 -case: H1=> t. 88 +by apply: or_introl. 89 +by apply: or_intror; apply: or_introl. 90 -by apply: or_intror; apply: or_intror. 91 -by apply: or_introl; apply: or_introl. 92 -case: H2=> t. 93 +by apply: or_introl; apply: or_intror. 94 +by apply: or_intror. 95 Qed Lemma myunioncompmother (A : myset M) : A (A^c) = mymotherset. 98 Proof. 99 apply: axiom_exteqmyset; rewrite / eqmyset / mysub; apply: conj => [x x HM] by case by case: ( axiom_myset A x); [ apply: or_introl apply: or_intror ]. 102 Qed. 103 End. mycupa myunioncompmother or_intror or_introl Definition mymap {M1 M2 : Type} (A : myset M1) (B : myset M2) 106 (f : M1 -> M2) 107 := (forall (x : M1), (x A) -> ((f x) B)). 108 Notation "f Map A \to B" := (mymap A B f) (at level 11).

29 'H 204 Abort 113 About 104 addn 43 addn1 44 addnc 45 Admitted 114 and 57, 76 apply/ 89 apply: 36, 73 apply: => 73 apply=> 73 Axiom 116 by 32 Canonical 120 case 58 case: 60 case => 59 case/ 90 case=> [ ] 78 Check 37, 103 CoInductive 201 Compute 102 coqc 204 Corollary 101 Defined 101 Definition 100 do 201 elim 79 End 32, 64 eq 43 exists 77, 123 Fact 101 field 201 Fixpoint 47, 101 Goal 56 H2 204 have 98 Hypothesis 29, 115 if 47 implicit 46 Inductive 42, 117 left 123 Lemma 101 Locate 110 Ltac 201 match with 43 move=> // 48 move/ 87 move: 31, 70 move: => 71 move=> 36, 69 move/ 55 Nat.add 43 O 42 or 76 Print 42, 105 Proof 31, 101 Proposition 101 Qed 32, 101 R 200 Record 118 Remark 101 Require Import 28, 205 rewrite 44, 82 rewrite /= 83 rewrite ( : = ) 49 rewrite / 54 right 123 S 42 Search 105 Section 28 Shift Ctrl C 44 Shift Ctrl P 41 split 123 suff 98 sum 47 Theorem 30, 101 Variable 114 wlog: 99 bigop 150 eqtype 131 fingroup 184, 192 finset 169 fintype 146, 166 Infotheo 196 Reals 200 seq 138 ssrbool 76, 126 ssrfun 46 ssrnat 41, 134 bool 75, 92 eqtype 131 False 77 list 124 nat 41, 77 Prop 29, 92, 117 seq 138 Set 117, 174 True 77 Type 117.vo AUTOMATH 10 Calculus of Constructions 14 Calculus of Inductive Constructions 14 CompCert 23 Coq 2 Coq/SSReflect/MathComp 2

30 211 CoqIDE 23 Coq 23 Display Notations 42 emacs 23 Gallina 14 itext4capofchans 203 MathComp 4 modus ponens 10 Open Scope 184 SSReflect 2 subgoal 30 System F , , , 42, 74, , 3, , 30 26, , , , , , 31, , 7 2, , , , ,

31 /4 2012/3 Research Scholar 2011/3 2012/ Reynald Affeldt 1976 = = 2000 Ingénieur Civil des Mines Coq/SSReflect/MathComp c FAX Printed in Japan ISBN

「計算と論理」 Software Foundations その4

「計算と論理」  Software Foundations   その4 Software Foundations 4 cal17@fos.kuis.kyoto-u.ac.jp http://www.fos.kuis.kyoto-u.ac.jp/~igarashi/class/cal/ November 7, 2017 ( ) ( 4) November 7, 2017 1 / 51 Poly.v ( ) ( 4) November 7, 2017 2 / 51 : (

More information

「計算と論理」 Software Foundations その3

「計算と論理」  Software Foundations   その3 Software Foundations 3 cal17@fos.kuis.kyoto-u.ac.jp October 24, 2017 ( ) ( 3) October 24, 2017 1 / 47 Lists.v ( ) ( ) ( ) ( 3) October 24, 2017 2 / 47 ( ) Inductive natprod : Type := pair : nat nat natprod.

More information

topics KNOPPIX/Math DVD maxima KSEG GeoGebra Coq 2011 July 17 - Page 1

topics KNOPPIX/Math DVD maxima KSEG GeoGebra Coq 2011 July 17 - Page 1 KNOPPIX/Math ( ) 2011/07/17 topics KNOPPIX/Math DVD maxima KSEG GeoGebra Coq 2011 July 17 - Page 1 (1) 2011 July 17 - Page 2 (2) 2011 July 17 - Page 3 KNOPPIX/Math KNOPPIX: Linux CD/DVD CD/DVD 1 Windows

More information

: Coq/SSReflect/MathComp, Coq., Coq SSReflect., MathComp,. Coq ( ) SSReflect, MathComp ( + ) :, Coq/SSReflect MathComp, : 1. Coq/SSReflect / / ( ) 2.

: Coq/SSReflect/MathComp, Coq., Coq SSReflect., MathComp,. Coq ( ) SSReflect, MathComp ( + ) :, Coq/SSReflect MathComp, : 1. Coq/SSReflect / / ( ) 2. @ 2015/7/24 2015 7 21( ) 24 ( ) : Coq/SSReflect/MathComp, Coq., Coq SSReflect., MathComp,. Coq ( ) SSReflect, MathComp ( + ) :, Coq/SSReflect MathComp, : 1. Coq/SSReflect / / ( ) 2. ( Coq ) 3. Coq SSReflect

More information

ML Edinburgh LCF ML Curry-Howard ML ( ) ( ) ( ) ( ) 1

ML Edinburgh LCF ML Curry-Howard ML ( ) ( ) ( ) ( ) 1 More Logic More Types ML/OCaml GADT Jacques Garrigue ( ) Jacques Le Normand (Google) Didier Rémy (INRIA) @garriguejej ocamlgadt ML Edinburgh LCF ML Curry-Howard ML ( ) ( ) ( ) ( ) 1 ( ) ML type nebou and

More information

Excel ではじめる数値解析 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

Excel ではじめる数値解析 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 初版 1 刷発行時のものです. Excel ではじめる数値解析 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/009631 このサンプルページの内容は, 初版 1 刷発行時のものです. Excel URL http://www.morikita.co.jp/books/mid/009631 i Microsoft Windows

More information

医系の統計入門第 2 版 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 第 2 版 1 刷発行時のものです.

医系の統計入門第 2 版 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 第 2 版 1 刷発行時のものです. 医系の統計入門第 2 版 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/009192 このサンプルページの内容は, 第 2 版 1 刷発行時のものです. i 2 t 1. 2. 3 2 3. 6 4. 7 5. n 2 ν 6. 2 7. 2003 ii 2 2013 10 iii 1987

More information

Akito Tsuboi June 22, T ϕ T M M ϕ M M ϕ T ϕ 2 Definition 1 X, Y, Z,... 1

Akito Tsuboi June 22, T ϕ T M M ϕ M M ϕ T ϕ 2 Definition 1 X, Y, Z,... 1 Akito Tsuboi June 22, 2006 1 T ϕ T M M ϕ M M ϕ T ϕ 2 Definition 1 X, Y, Z,... 1 1. X, Y, Z,... 2. A, B (A), (A) (B), (A) (B), (A) (B) Exercise 2 1. (X) (Y ) 2. ((X) (Y )) (Z) 3. (((X) (Y )) (Z)) Exercise

More information

<4D F736F F D B B BB2D834A836F815B82D082C88C602E646F63>

<4D F736F F D B B BB2D834A836F815B82D082C88C602E646F63> 入門モーター工学 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/074351 このサンプルページの内容は, 初版 1 刷発行当時のものです. 10 kw 21 20 50 2 20 IGBT IGBT IGBT 21 (1) 1 2 (2) (3) ii 20 2013 2 iii iv...

More information

koba/class/soft-kiso/ 1 λ if λx.λy.y false 0 λ typed λ-calculus λ λ 1.1 λ λ, syntax τ (types) ::= b τ 1 τ 2 τ 1

koba/class/soft-kiso/ 1 λ if λx.λy.y false 0 λ typed λ-calculus λ λ 1.1 λ λ, syntax τ (types) ::= b τ 1 τ 2 τ 1 http://www.kb.ecei.tohoku.ac.jp/ koba/class/soft-kiso/ 1 λ if λx.λy.y false 0 λ typed λ-calculus λ λ 1.1 λ 1.1.1 λ, syntax τ (types) ::= b τ 1 τ 2 τ 1 τ 2 M (terms) ::= c τ x M 1 M 2 λx : τ.m (M 1,M 2

More information

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63>

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63> デザイン言語 Processing 入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/084931 このサンプルページの内容は, 初版 1 刷発行当時のものです. Processing Ben Fry Casey Reas Windows Mac Linux Lesson 1 Processing

More information

<4D F736F F D B B BB2D834A836F815B82D082C88C60202D B2E646F63>

<4D F736F F D B B BB2D834A836F815B82D082C88C60202D B2E646F63> 例題で学ぶはじめての塑性力学 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/066721 このサンプルページの内容は, 初版 1 刷発行当時のものです. http://www.morikita.co.jp/support/ 03 3817 5670 FAX 03 3815 8199 i 1

More information

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63>

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63> 新 Excel コンピュータシミュレーション サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/084871 このサンプルページの内容は, 初版 1 刷発行当時のものです. Microsoft Excel Excel Visual Basic Visual Basic 2007 Excel Excel

More information

Objective Caml 3.12 Jacques Garrigue ( ) with Alain Frisch (Lexifi), OCaml developper team (INRIA)

Objective Caml 3.12 Jacques Garrigue ( )   with Alain Frisch (Lexifi), OCaml developper team (INRIA) Objective Caml 3.12 Jacques Garrigue ( ) http://www.math.nagoya-u.ac.jp/~garrigue/ with Alain Frisch (Lexifi), OCaml developper team (INRIA) Jacques Garrigue Modules in Objective Caml 3.12 1 Objective

More information

Copyright c 2008 Zhenjiang Hu, All Right Reserved.

Copyright c 2008 Zhenjiang Hu, All Right Reserved. 2008 10 27 Copyright c 2008 Zhenjiang Hu, All Right Reserved. (Bool) True False data Bool = False True Remark: not :: Bool Bool not False = True not True = False (Pattern matching) (Rewriting rules) not

More information

微分積分 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

微分積分 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 初版 1 刷発行時のものです. 微分積分 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. ttp://www.morikita.co.jp/books/mid/00571 このサンプルページの内容は, 初版 1 刷発行時のものです. i ii 014 10 iii [note] 1 3 iv 4 5 3 6 4 x 0 sin x x 1 5 6 z = f(x, y) 1 y = f(x)

More information

newmain.dvi

newmain.dvi 数論 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/008142 このサンプルページの内容は, 第 2 版 1 刷発行当時のものです. Daniel DUVERNEY: THÉORIE DES NOMBRES c Dunod, Paris, 1998, This book is published

More information

I: 2 : 3 +

I: 2 : 3 + I: 1 I: 2008 I: 2 : 3 + I: 3, 3700. (ISBN4-00-010352-0) H.P.Barendregt, The lambda calculus: its syntax and semantics, Studies in logic and the foundations of mathematics, v.103, North-Holland, 1984. (ISBN

More information

provider_020524_2.PDF

provider_020524_2.PDF 1 1 1 2 2 3 (1) 3 (2) 4 (3) 6 7 7 (1) 8 (2) 21 26 27 27 27 28 31 32 32 36 1 1 2 2 (1) 3 3 4 45 (2) 6 7 5 (3) 6 7 8 (1) ii iii iv 8 * 9 10 11 9 12 10 13 14 15 11 16 17 12 13 18 19 20 (2) 14 21 22 23 24

More information

Parametric Polymorphism

Parametric Polymorphism ML 2 2011/04/19 Parametric Polymorphism Type Polymorphism ? : val hd_int : int list - > int val hd_bool : bool list - > bool val hd_i_x_b : (int * bool) list - > int * bool etc. let hd_int = function (x

More information

44 4 I (1) ( ) (10 15 ) ( 17 ) ( 3 1 ) (2)

44 4 I (1) ( ) (10 15 ) ( 17 ) ( 3 1 ) (2) (1) I 44 II 45 III 47 IV 52 44 4 I (1) ( ) 1945 8 9 (10 15 ) ( 17 ) ( 3 1 ) (2) 45 II 1 (3) 511 ( 451 1 ) ( ) 365 1 2 512 1 2 365 1 2 363 2 ( ) 3 ( ) ( 451 2 ( 314 1 ) ( 339 1 4 ) 337 2 3 ) 363 (4) 46

More information

i ii i iii iv 1 3 3 10 14 17 17 18 22 23 28 29 31 36 37 39 40 43 48 59 70 75 75 77 90 95 102 107 109 110 118 125 128 130 132 134 48 43 43 51 52 61 61 64 62 124 70 58 3 10 17 29 78 82 85 102 95 109 iii

More information

# let st1 = {name = "Taro Yamada"; id = };; val st1 : student = {name="taro Yamada"; id=123456} { 1 = 1 ;...; n = n } # let string_of_student {n

# let st1 = {name = Taro Yamada; id = };; val st1 : student = {name=taro Yamada; id=123456} { 1 = 1 ;...; n = n } # let string_of_student {n II 6 / : 2001 11 21 (OCaml ) 1 (field) name id type # type student = {name : string; id : int};; type student = { name : string; id : int; } student {} type = { 1 : 1 ;...; n : n } { 1 = 1 ;...; n = n

More information

Copyright c 2006 Zhenjiang Hu, All Right Reserved.

Copyright c 2006 Zhenjiang Hu, All Right Reserved. 1 2006 Copyright c 2006 Zhenjiang Hu, All Right Reserved. 2 ( ) 3 (T 1, T 2 ) T 1 T 2 (17.3, 3) :: (Float, Int) (3, 6) :: (Int, Int) (True, (+)) :: (Bool, Int Int Int) 4 (, ) (, ) :: a b (a, b) (,) x y

More information

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C602E646F63>

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C602E646F63> スピントロニクスの基礎 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/077461 このサンプルページの内容は, 初版 1 刷発行時のものです. i 1 2 ii 3 5 4 AMR (anisotropic magnetoresistance effect) GMR (giant magnetoresistance

More information

# let rec sigma (f, n) = # if n = 0 then 0 else f n + sigma (f, n-1);; val sigma : (int -> int) * int -> int = <fun> sigma f n ( : * -> * ) sqsum cbsu

# let rec sigma (f, n) = # if n = 0 then 0 else f n + sigma (f, n-1);; val sigma : (int -> int) * int -> int = <fun> sigma f n ( : * -> * ) sqsum cbsu II 4 : 2001 11 7 keywords: 1 OCaml OCaml (first-class value) (higher-order function) 1.1 1 2 + 2 2 + + n 2 sqsum 1 3 + 2 3 + + n 3 cbsum # let rec sqsum n = # if n = 0 then 0 else n * n + sqsum (n - 1)

More information

; Modus Ponens 1

; Modus Ponens 1 1 9 00 ; 1402 5 16 20 1502 1 11 1 1 2 1 2 Modus Ponens 1 1 2 Modus Ponens 2 1 12 Gentzen 13 Modus ponens 1 100 2 100 100 P Q P Q Q 2 P Q P Q Modus ponens Y Y 1 Modus Ponens P 2 Y Y Y Y Y Y C D Y F (C D)

More information

地盤環境振動の対策技術-00-前付.indd

地盤環境振動の対策技術-00-前付.indd 地盤環境振動の対策技術 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/048561 このサンプルページの内容は, 初版 1 刷発行当時のものです. i 23 25 28 8 ii 1 8 2 9 3 10 4 11 5 12 6 13 7 iii 1 1 1.1 1.1.11 1.1.22

More information

Jacques Garrigue

Jacques Garrigue Jacques Garrigue Garrigue 1 Garrigue 2 $ print_lines () > for i in $1; do > echo $i > done $ print_lines "a b c" a b c Garrigue 3 Emacs Lisp (defun print-lines (lines) (dolist (str lines) (insert str)

More information

論理学入門 講義ノート email: mitsu@abelardfletkeioacjp Copyright c 1995 by the author ll right reserved 1 1 3 2 5 3 7 31 7 32 9 33 13 4 29 41 33 42 38 5 45 51 45 52 47 3 1 19 [ 1] Begin at the beginning [ 2] [

More information

JavaCard p.1/41

JavaCard   p.1/41 JavaCard Email : nagamiya@comp.cs.gunma-u.ac.jp p.1/41 Hoare Java p.2/41 (formal method) (formal specification) (formal) JML, D, VDM, (formal method) p.3/41 Hoare Java p.4/41 (precondition) (postcondition)

More information

フリーソフトでつくる音声認識システム ( 第 2 版 ) サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 第 2 版 1 刷発行時のものです.

フリーソフトでつくる音声認識システム ( 第 2 版 ) サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 第 2 版 1 刷発行時のものです. フリーソフトでつくる音声認識システム ( 第 2 版 ) サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/084712 このサンプルページの内容は, 第 2 版 1 刷発行時のものです. i 2007 10 1 Scilab 2 2017 2 1 2 1 ii 2 web 2007 9 iii

More information

数理計画法入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

数理計画法入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 初版 1 刷発行時のものです. 数理計画法入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/092181 このサンプルページの内容は, 初版 1 刷発行時のものです. i 1947 G.B. Dantzig 3 (1) (2) (3) (4) Microsoft Excel Web 4 1 2 2 2 2 3 ii 4

More information

例題で学ぶオペレーションズ リサーチ入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

例題で学ぶオペレーションズ リサーチ入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 初版 1 刷発行時のものです. 例題で学ぶオペレーションズ リサーチ入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/009641 このサンプルページの内容は, 初版 1 刷発行時のものです. i OR OR OR OR OR OR OR OR OR 2015 5 ii 1 OR 1 1.1 OR... 1 1.2 OR...

More information

VDM-SL VDM VDM-SL Toolbox VDM++ Toolbox 1 VDM-SL VDM++ Web bool

VDM-SL VDM VDM-SL Toolbox VDM++ Toolbox 1 VDM-SL VDM++ Web bool VDM-SL VDM++ 23 6 28 VDM-SL Toolbox VDM++ Toolbox 1 VDM-SL VDM++ Web 2 1 3 1.1............................................... 3 1.1.1 bool......................................... 3 1.1.2 real rat int

More information

SCM (v0201) ( ) SCM 2 SCM 3 SCM SCM 2.1 SCM SCM SCM (1) MS-DOS (2) Microsoft(R) Windows 95 (C)Copyright Microsoft Corp

SCM (v0201) ( ) SCM 2 SCM 3 SCM SCM 2.1 SCM SCM SCM (1) MS-DOS (2) Microsoft(R) Windows 95 (C)Copyright Microsoft Corp SCM (v0201) ( ) 14 4 20 1 SCM 2 SCM 3 SCM 4 5 2 SCM 2.1 SCM SCM 2 1 2 SCM (1) MS-DOS (2) Microsoft(R) Windows 95 (C)Copyright Microsoft Corp 1981-1996. 1 (3) C:\WINDOWS>cd.. C:\>cd scm C:\SCM> C:\SCM>

More information

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63>

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63> 常微分方程式の局所漸近解析 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/007651 このサンプルページの内容は, 初版 1 刷発行当時のものです. i Leibniz ydy = y 2 /2 1675 11 11 [6] 100 Bernoulli Riccati 19 Fuchs

More information

並列計算の数理とアルゴリズム サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

並列計算の数理とアルゴリズム サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.  このサンプルページの内容は, 初版 1 刷発行時のものです. 並列計算の数理とアルゴリズム サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/080711 このサンプルページの内容は, 初版 1 刷発行時のものです. Calcul scientifique parallèle by Frédéric Magoulès and François-Xavier

More information

Int Int 29 print Int fmt tostring 2 2 [19] ML ML [19] ML Emacs Standard ML M M ::= x c λx.m M M let x = M in M end (M) x c λx.

Int Int 29 print Int fmt tostring 2 2 [19] ML ML [19] ML Emacs Standard ML M M ::= x c λx.m M M let x = M in M end (M) x c λx. 1, 2 1 m110057@shibaura-it.ac.jp 2 sasano@sic.shibaura-it.ac.jp Eclipse Visual Studio ML Standard ML Emacs 1 ( IDE ) IDE C C++ Java IDE IDE IDE IDE Eclipse Java IDE Java Standard ML 1 print (Int. 1 Int

More information

25 II :30 16:00 (1),. Do not open this problem booklet until the start of the examination is announced. (2) 3.. Answer the following 3 proble

25 II :30 16:00 (1),. Do not open this problem booklet until the start of the examination is announced. (2) 3.. Answer the following 3 proble 25 II 25 2 6 13:30 16:00 (1),. Do not open this problem boolet until the start of the examination is announced. (2) 3.. Answer the following 3 problems. Use the designated answer sheet for each problem.

More information

Tricorn

Tricorn Triorn 016 3 1 Mandelbrot Triorn Mandelbrot Robert L DevaneyAn introdution to haoti dynamial Systems Addison-Wesley, 1989 Triorn 1 W.D.Crowe, R.Hasson, P.J.Rippon, P.E.D.Strain- Clark, On the struture

More information

org/ghc/ Windows Linux RPM 3.2 GHCi GHC gcc javac ghc GHCi(ghci) GHCi Prelude> GHCi :load file :l file :also file :a file :reload :r :type expr :t exp

org/ghc/ Windows Linux RPM 3.2 GHCi GHC gcc javac ghc GHCi(ghci) GHCi Prelude> GHCi :load file :l file :also file :a file :reload :r :type expr :t exp 3 Haskell Haskell Haskell 1. 2. 3. 4. 5. 1. 2. 3. 4. 5. 6. C Java 3.1 Haskell Haskell GHC (Glasgow Haskell Compiler 1 ) GHC Haskell GHC http://www.haskell. 1 Guarded Horn Clauses III - 1 org/ghc/ Windows

More information

untitled

untitled Trademark of American Soybean Association TM http://www.wakachiku.co.jp 8080024 147 TEL 0937611331 1530064 22318 TEL 0334920271 0640807 1136 2 TEL 0115111881 9800014 21028 TEL 0222214325 2600022 322 TEL

More information

MS55D_J

MS55D_J POWERED MULTIMEDIA SPEAKERS 0 10 YST-MS55D POWERED MULTIMEDIA SPEAKERS VOLUME YST-MS55D POWERED MULTIMEDIA SPEAKERS BASS ii iii iv POWERED MULTIMEDIA SPEAKERS YST-MS55D BASS 0 10 POWERED MULTIMEDIA SPEAKERS

More information

Test IV, March 22, 2016 6. Suppose that 2 n a n converges. Prove or disprove that a n converges. Proof. Method I: Let a n x n be a power series, which converges at x = 2 by the assumption. Applying Theorem

More information

ルベーグ積分 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 初版 1 刷発行時のものです.

ルベーグ積分 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.   このサンプルページの内容は, 初版 1 刷発行時のものです. ルベーグ積分 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/005431 このサンプルページの内容は, 初版 1 刷発行時のものです. Lebesgue 1 2 4 4 1 2 5 6 λ a

More information

Emacs Ruby..

Emacs Ruby.. command line editor 27014533 2018 3 1 5 1.1................................... 5 1.2................................... 5 2 6 2.1 Emacs...................................... 6 2.2 Ruby.......................................

More information

haskell.gby

haskell.gby Haskell 1 2 3 Haskell ( ) 4 Haskell Lisper 5 Haskell = Haskell 6 Haskell Haskell... 7 qsort [8,2,5,1] [1,2,5,8] "Hello, " ++ "world!" "Hello, world!" 1 + 2 div 8 2 (+) 1 2 8 div 2 3 4 map even [1,2,3,4]

More information

=

= 2. 2.1 2.2 kuri@ice.uec.ac.jp ( 2007/10/30/16:46) 1 . 1. 1 + 2 = 5. 2. 180. 3. 3 3. 4.. 5.. 2 2.1 1.,,,,. 2., ( ) ( ).,,,, 3.,. 4.,,,. 3 1.,. 1. 1 + 2 = 5. (, ) 2. 180. (, ) 3. 3, 3. (, ) 4.. (, ) 5..

More information

2

2 01 02 03 04 05 06 07 08 09 10 11 12 13 14 15 16 17 18 19 20 21 22 23 24 2 3 01 02 03 4 04 05 06 5 07 08 09 6 10 11 12 7 13 14 15 8 16 17 18 9 19 20 21 10 22 23 24 11 FIELD MAP 12 13 http://www.pref.ishikawa.jp/shinrin/zei/index.html

More information

0.2 Button TextBox: menu tab 2

0.2 Button TextBox: menu tab 2 Specview VO 2012 2012/9/27 Specview Specview STSCI(Space Telescope SCience Institute) VO Specview Web page http://www.stsci.edu/resources/software hardware/specview http://specview.stsci.edu/javahelp/main.html

More information

i

i 14 i ii iii iv v vi 14 13 86 13 12 28 14 16 14 15 31 (1) 13 12 28 20 (2) (3) 2 (4) (5) 14 14 50 48 3 11 11 22 14 15 10 14 20 21 20 (1) 14 (2) 14 4 (3) (4) (5) 12 12 (6) 14 15 5 6 7 8 9 10 7

More information

( ) P, P P, P (negation, NOT) P ( ) P, Q, P Q, P Q 3, P Q (logical product, AND) P Q ( ) P, Q, P Q, P Q, P Q (logical sum, OR) P Q ( ) P, Q, P Q, ( P

( ) P, P P, P (negation, NOT) P ( ) P, Q, P Q, P Q 3, P Q (logical product, AND) P Q ( ) P, Q, P Q, P Q, P Q (logical sum, OR) P Q ( ) P, Q, P Q, ( P Advent Calendar 2018 @Fukuso Sutaro,,, ( ) Davidson, 5, 1 (quantification) (open sentence) 1,,,,,, 1 1 (propositional logic) (truth value) (proposition) (sentence) 2 (2-valued logic) 2, true false (truth

More information

II

II II 2016 7 21 computer-assisted proof 1 / 64 1. 2. 3. Siegfried M. Rump : [1] I,, 14:3 (2004), pp. 214 223. [2] II,, 14:4 (2004), pp. 346 359. 2 / 64 Risch 18 3 / 64 M n = 2 n 1 (n = 1, 2,... ) 2 2 1 1

More information

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63>

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63> 電気電子数学入門 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/073471 このサンプルページの内容は, 初版 1 刷発行当時のものです. i 14 (tool) [ ] IT ( ) PC (EXCEL) HP() 1 1 4 15 3 010 9 ii 1... 1 1.1 1 1.

More information

( ) ( ) lex LL(1) LL(1)

( ) ( ) lex LL(1) LL(1) () () lex LL(1) LL(1) http://www.cs.info.mie-u.ac.jp/~toshi/lectures/compiler/ 29 5 14 1 1 () / (front end) (back end) (phase) (pass) 1 2 1 () () var left, right; fun int main() { left = 0; right = 10;

More information

fp.gby

fp.gby 1 1 2 2 3 2 4 5 6 7 8 9 10 11 Haskell 12 13 Haskell 14 15 ( ) 16 ) 30 17 static 18 (IORef) 19 20 OK NG 21 Haskell (+) :: Num a => a -> a -> a sort :: Ord a => [a] -> [a] delete :: Eq a => a -> [a] -> [a]

More information

第1部 一般的コメント

第1部 一般的コメント (( 2000 11 24 2003 12 31 3122 94 2332 508 26 a () () i ii iii iv (i) (ii) (i) (ii) (iii) (iv) (a) (b)(c)(d) a) / (i) (ii) (iii) (iv) 1996 7 1996 12

More information

表1票4.qx4

表1票4.qx4 iii iv v 2 3 4 5 6 7 8 9 10 11 12 13 14 15 16 17 18 19 22 23 10 11 24 25 26 27 10 56 28 11 29 30 12 13 14 15 16 17 18 19 2010 2111 22 23 2412 2513 14 31 17 32 18 33 19 34 20 35 21 36 24 37 25 38 2614

More information

HARK Designer Documentation 0.5.0 HARK support team 2013 08 13 Contents 1 3 2 5 2.1.......................................... 5 2.2.............................................. 5 2.3 1: HARK Designer.................................

More information

第1章 国民年金における無年金

第1章 国民年金における無年金 1 2 3 4 ILO ILO 5 i ii 6 7 8 9 10 ( ) 3 2 ( ) 3 2 2 2 11 20 60 12 1 2 3 4 5 6 7 8 9 10 11 12 13 13 14 15 16 17 14 15 8 16 2003 1 17 18 iii 19 iv 20 21 22 23 24 25 ,,, 26 27 28 29 30 (1) (2) (3) 31 1 20

More information

C による数値計算法入門 ( 第 2 版 ) 新装版 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. このサンプルページの内容は, 新装版 1 刷発行時のものです.

C による数値計算法入門 ( 第 2 版 ) 新装版 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます.  このサンプルページの内容は, 新装版 1 刷発行時のものです. C による数値計算法入門 ( 第 2 版 ) 新装版 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/009383 このサンプルページの内容は, 新装版 1 刷発行時のものです. i 2 22 2 13 ( ) 2 (1) ANSI (2) 2 (3) Web http://www.morikita.co.jp/books/mid/009383

More information

GNU Emacs GNU Emacs

GNU Emacs GNU Emacs GNU Emacs 2015 10 2 1 GNU Emacs 1 1.1....................................... 1 1.2....................................... 1 1.2.1..................................... 1 1.2.2.....................................

More information

New version (2.15.1) of Specview is now available Dismiss Windows Specview.bat set spv= Specview set jhome= JAVA (C:\Program Files\Java\jre<version>\

New version (2.15.1) of Specview is now available Dismiss Windows Specview.bat set spv= Specview set jhome= JAVA (C:\Program Files\Java\jre<version>\ Specview VO 2012 2012/3/26 Specview Specview STSCI(Space Telescope SCience Institute) VO Specview Web page http://www.stsci.edu/resources/software hardware/specview http://specview.stsci.edu/javahelp/main.html

More information

コンピュータ概論

コンピュータ概論 4.1 For Check Point 1. For 2. 4.1.1 For (For) For = To Step (Next) 4.1.1 Next 4.1.1 4.1.2 1 i 10 For Next Cells(i,1) Cells(1, 1) Cells(2, 1) Cells(10, 1) 4.1.2 50 1. 2 1 10 3. 0 360 10 sin() 4.1.2 For

More information

<4D F736F F D B B BB2D834A836F815B82D082C88C602E646F63>

<4D F736F F D B B BB2D834A836F815B82D082C88C602E646F63> 信号処理の基礎 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/081051 このサンプルページの内容は, 初版 1 刷発行時のものです. i AI ii z / 2 3 4 5 6 7 7 z 8 8 iii 2013 3 iv 1 1 1.1... 1 1.2... 2 2 4 2.1...

More information

X Window System X X &

X Window System X X & 1 1 1.1 X Window System................................... 1 1.2 X......................................... 1 1.3 X &................................ 1 1.3.1 X.......................... 1 1.3.2 &....................................

More information

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63>

<4D F736F F D B B83578B6594BB2D834A836F815B82D082C88C60202E646F63> 単純適応制御 SAC サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/091961 このサンプルページの内容は, 初版 1 刷発行当時のものです. 1 2 3 4 5 9 10 12 14 15 A B F 6 8 11 13 E 7 C D URL http://www.morikita.co.jp/support

More information

<4D F736F F D B B BB2D834A836F815B82D082C88C60202D B2E646F63>

<4D F736F F D B B BB2D834A836F815B82D082C88C60202D B2E646F63> 入社 5 年目までに身につけたい建設エンジニアの仕事術 サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/087141 このサンプルページの内容は, 初版 1 刷発行当時のものです. i 3 5 2009 1 ii 1 1 1 2 3 3 6 13 1.1 14 1.2 15 1.3 17 1.4

More information

20 15 14.6 15.3 14.9 15.7 16.0 15.7 13.4 14.5 13.7 14.2 10 10 13 16 19 22 1 70,000 60,000 50,000 40,000 30,000 20,000 10,000 0 2,500 59,862 56,384 2,000 42,662 44,211 40,639 37,323 1,500 33,408 34,472

More information

- 2 -

- 2 - - 2 - - 3 - (1) (2) (3) (1) - 4 - ~ - 5 - (2) - 6 - (1) (1) - 7 - - 8 - (i) (ii) (iii) (ii) (iii) (ii) 10 - 9 - (3) - 10 - (3) - 11 - - 12 - (1) - 13 - - 14 - (2) - 15 - - 16 - (3) - 17 - - 18 - (4) -

More information

2 1980 8 4 4 4 4 4 3 4 2 4 4 2 4 6 0 0 6 4 2 4 1 2 2 1 4 4 4 2 3 3 3 4 3 4 4 4 4 2 5 5 2 4 4 4 0 3 3 0 9 10 10 9 1 1

2 1980 8 4 4 4 4 4 3 4 2 4 4 2 4 6 0 0 6 4 2 4 1 2 2 1 4 4 4 2 3 3 3 4 3 4 4 4 4 2 5 5 2 4 4 4 0 3 3 0 9 10 10 9 1 1 1 1979 6 24 3 4 4 4 4 3 4 4 2 3 4 4 6 0 0 6 2 4 4 4 3 0 0 3 3 3 4 3 2 4 3? 4 3 4 3 4 4 4 4 3 3 4 4 4 4 2 1 1 2 15 4 4 15 0 1 2 1980 8 4 4 4 4 4 3 4 2 4 4 2 4 6 0 0 6 4 2 4 1 2 2 1 4 4 4 2 3 3 3 4 3 4 4

More information

I? 3 1 3 1.1?................................. 3 1.2?............................... 3 1.3!................................... 3 2 4 2.1........................................ 4 2.2.......................................

More information

1 (1) (2)

1 (1) (2) 1 2 (1) (2) (3) 3-78 - 1 (1) (2) - 79 - i) ii) iii) (3) (4) (5) (6) - 80 - (7) (8) (9) (10) 2 (1) (2) (3) (4) i) - 81 - ii) (a) (b) 3 (1) (2) - 82 - - 83 - - 84 - - 85 - - 86 - (1) (2) (3) (4) (5) (6)

More information

main.dvi

main.dvi Java でつくる RoboCup サッカー選手プログラム サンプルページ この本の定価 判型などは, 以下の URL からご覧いただけます. http://www.morikita.co.jp/books/mid/084531 このサンプルページの内容は, 初版 1 刷発行当時のものです. http://www.morikita.co.jp/soft/robocup/ ( 03 3817 5670

More information

T rank A max{rank Q[R Q, J] t-rank T [R T, C \ J] J C} 2 ([1, p.138, Theorem 4.2.5]) A = ( ) Q rank A = min{ρ(j) γ(j) J J C} C, (5) ρ(j) = rank Q[R Q,

T rank A max{rank Q[R Q, J] t-rank T [R T, C \ J] J C} 2 ([1, p.138, Theorem 4.2.5]) A = ( ) Q rank A = min{ρ(j) γ(j) J J C} C, (5) ρ(j) = rank Q[R Q, (ver. 4:. 2005-07-27) 1 1.1 (mixed matrix) (layered mixed matrix, LM-matrix) m n A = Q T (2m) (m n) ( ) ( ) Q I m Q à = = (1) T diag [t 1,, t m ] T rank à = m rank A (2) 1.2 [ ] B rank [B C] rank B rank

More information

18 5 10 1 1 1.1 1.1.1 P Q P Q, P, Q P Q P Q P Q, P, Q 2 1 1.1.2 P.Q T F Z R 0 1 x, y x + y x y x y = y x x (y z) = (x y) z x + y = y + x x + (y + z) = (x + y) + z P.Q V = {T, F } V P.Q P.Q T F T F 1.1.3

More information

Excel97関数編

Excel97関数編 Excel97 SUM Microsoft Excel 97... 1... 1... 1... 2... 3... 3... 4... 5... 6... 6... 7 SUM... 8... 11 Microsoft Excel 97 AVERAGE MIN MAX SUM IF 2 RANK TODAY ROUND COUNT INT VLOOKUP 1/15 Excel A B C A B

More information

Introduction Purpose This training course demonstrates the use of the High-performance Embedded Workshop (HEW), a key tool for developing software for

Introduction Purpose This training course demonstrates the use of the High-performance Embedded Workshop (HEW), a key tool for developing software for Introduction Purpose This training course demonstrates the use of the High-performance Embedded Workshop (HEW), a key tool for developing software for embedded systems that use microcontrollers (MCUs)

More information

III III 2010 PART I 1 Definition 1.1 (, σ-),,,, Borel( ),, (σ-) (M, F, µ), (R, B(R)), (C, B(C)) Borel Definition 1.2 (µ-a.e.), (in µ), (in L 1 (µ)). T

III III 2010 PART I 1 Definition 1.1 (, σ-),,,, Borel( ),, (σ-) (M, F, µ), (R, B(R)), (C, B(C)) Borel Definition 1.2 (µ-a.e.), (in µ), (in L 1 (µ)). T III III 2010 PART I 1 Definition 1.1 (, σ-),,,, Borel( ),, (σ-) (M, F, µ), (R, B(R)), (C, B(C)) Borel Definition 1.2 (µ-a.e.), (in µ), (in L 1 (µ)). Theorem 1.3 (Lebesgue ) lim n f n = f µ-a.e. g L 1 (µ)

More information

Microsoft PowerPoint - ProD0107.ppt

Microsoft PowerPoint - ProD0107.ppt プログラミング D M 講義資料 教科書 :6 章 中田明夫 nakata@ist.osaka-u.ac.jp 2005/1/7 プログラミング D -M- 1 2005/1/7 プログラミング D -M- 2 リスト 1 リスト : 同じ型の値の並び val h=[10,6,7,8,~8,5,9]; val h = [10,6,7,8,~8,5,9]: int list val g=[1.0,4.5,

More information

パズルをSugar制約ソルバーで解く

パズルをSugar制約ソルバーで解く Sugar 1 2 3 1 CSPSAT 2008 8 21 Sugar 1 2 3 Sugar Sugar (CSP) (SAT ) (encode) SAT SAT order encoding direct encoding support encoding http://bachistckobe-uacjp/sugar/ Web Sugar 1 2 3 Sugar SAT (COP) MAX-CSP

More information

1st-session key

1st-session key 1 2013/11/29 Project based Learning: Soccer Agent Program 1 2012/12/9 Project based Learning: Soccer Agent Program PBL Learning by doing Schedule 1,2 2013 11/29 Make 2013 12/6 2013 12/13 2013 12/20 2014

More information

Specview Specview Specview STSCI(Space Telescope SCience Institute) VO Specview Web page htt

Specview Specview Specview STSCI(Space Telescope SCience Institute) VO Specview Web page   htt Specview Specview Specview STSCI(Space Telescope SCience Institute) VO Specview Web page http://www.stsci.edu/resources/software_hardware/specview http://specview.stsci.edu/javahelp/main.html Specview

More information

syspro-0405.ppt

syspro-0405.ppt 3 4, 5 1 UNIX csh 2.1 bash X Window 2 grep l POSIX * more POSIX 3 UNIX. 4 first.sh #!bin/sh #first.sh #This file looks through all the files in the current #directory for the string yamada, and then prints

More information

RQT8189-S.indd

RQT8189-S.indd A Operating Instructions Portable CD Player SL-CT730 BATTERY CARRYING CASE SL-CT730 SL-CT830 RQT8189-S F0805SZ0 OPEN OPEN + - + - DC IN SL-CT730SL-CT830 DC IN EXT BATT DC IN () SL-CT730 SL-CT830 SL-CT730

More information

橡最新卒論

橡最新卒論 Research of improving of recognition ability in Face recognition system Abstract The age when baiometrics was used as a password came today. Because various baiometrics such as a voice, a fingerprint,

More information